Skip to content

Commit

Permalink
chore: improve doc string
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Jan 9, 2025
1 parent de2f4e2 commit c5282db
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Grind/Offset.lean
Original file line number Diff line number Diff line change
Expand Up @@ -126,7 +126,7 @@ theorem Cnstrs.unsat' (ctx : Context) (c : Cnstrs) : c.isFalse = true → ¬ c.d
have := Cnstr.of_isFalse ctx h₁
contradiction

/-- Returns `c_1 → ... → c_n → C -/
/-- `denote ctx [c_1, ..., c_n] C` is `c_1.denote ctx → ... → c_n.denote ctx → C` -/
def Cnstrs.denote (ctx : Context) (cs : Cnstrs) (C : Prop) : Prop :=
match cs with
| [] => C
Expand Down

0 comments on commit c5282db

Please sign in to comment.