Skip to content

Commit

Permalink
checkpoint
Browse files Browse the repository at this point in the history
  • Loading branch information
markusdemedeiros committed Nov 5, 2024
1 parent 81ecab6 commit fd2fb82
Showing 1 changed file with 15 additions and 0 deletions.
15 changes: 15 additions & 0 deletions SampCert/Foundations/While.lean
Original file line number Diff line number Diff line change
Expand Up @@ -58,4 +58,19 @@ theorem probWhile_apply (cond : T → Bool) (body : T → SLang T) (init : T) (x
· apply probWhileCut_monotonic
· apply H


-- A version of probWhile that proves normalization, when its arguments are all normal
def SPMF_while (cond : T → Bool) (body : T → SPMF T) (init : T) : SPMF T :=
⟨ probWhile cond (fun x => body x) init,
by
unfold probWhile
sorry

lemma SPMF_while_eq (cond : T → Bool) (body : T → SPMF T) (init : T) :
((SPMF_while cond body init) : SLang T) = (probWhile cond (fun x => body x) init) := by
simp [SPMF_while]




end SLang

0 comments on commit fd2fb82

Please sign in to comment.