Skip to content

Commit

Permalink
start with "starCases"
Browse files Browse the repository at this point in the history
  • Loading branch information
m4lvin committed Oct 18, 2023
1 parent 07f9d0e commit d84f57e
Show file tree
Hide file tree
Showing 2 changed files with 17 additions and 1 deletion.
17 changes: 16 additions & 1 deletion Pdl/Semantics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,14 +22,29 @@ inductive StarCat {α : Type} (r : α → α → Prop) : α → α → Prop
| refl (a : α) : StarCat r a a
| step (a b c : α) : r a b → StarCat r b c → StarCat r a c


theorem StarIncl {α : Type} {a : α} {b : α} {r : α → α → Prop} : r a b → StarCat r a b :=
by
intro a_r_b
apply StarCat.step
exact a_r_b
exact StarCat.refl b

theorem starCases {α : Type} {a c : α} {r : α → α → Prop} :
StarCat r a c ↔ a = c ∨ (a ≠ c ∧ ∃ b, r a b ∧ StarCat r b c) :=
by
constructor
· intro r_aS_c
sorry
· intro rhs
cases rhs
case inl a_is_c =>
subst a_is_c
apply StarCat.refl
case inr hyp =>
rcases hyp with ⟨_, b, b_aS_c⟩
apply StarCat.step a b c
tauto
tauto
mutual
@[simp]
def evaluate {W : Type} : KripkeModel W → W → Formula → Prop
Expand Down
1 change: 1 addition & 0 deletions Pdl/Unravel.lean
Original file line number Diff line number Diff line change
Expand Up @@ -223,6 +223,7 @@ theorem likeLemmaFour :
absurd w_neq_v
rfl
case step u w_a_u u_aS_v =>
-- idea: use starCases here?
have IHa := likeLemmaFour M a w u X'
specialize IHa (⌈∗a⌉P) _ _ w_a_u _
· sorry
Expand Down

0 comments on commit d84f57e

Please sign in to comment.