Skip to content

Commit

Permalink
修正
Browse files Browse the repository at this point in the history
  • Loading branch information
Seasawher committed Oct 8, 2024
1 parent 67f4988 commit 3436d7f
Showing 1 changed file with 3 additions and 5 deletions.
8 changes: 3 additions & 5 deletions ConcreteSemantics/EquivalenceWithBigStep.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ BigStep 意味論を、SmallStep に翻訳できる。
-/
import ConcreteSemantics.BigStep
import ConcreteSemantics.SmallStep
import Mathlib.Tactic

open Relation

Expand All @@ -23,11 +22,10 @@ theorem big_step_to_small_step_star {S : Stmt} {s t : State} (h : (S, s) ==> t)
_ ⇒* (_, _) := by small_step

case step1 =>
set ct := (skip, t₁) with hcs
generalize hct : (skip, t₁) = ct
rw [hct] at hS_ih
induction hS_ih
case refl => rfl
case refl => sorry
case tail _ _ _ =>

sorry
-- apply SmallStep.seq_step (hS := hS₁)
sorry

0 comments on commit 3436d7f

Please sign in to comment.