Skip to content

Commit

Permalink
fix(data/fintype/basic): move card_subtype_mono into the fintype name…
Browse files Browse the repository at this point in the history
…space (#15185)
  • Loading branch information
linesthatinterlace committed Jul 8, 2022
1 parent 1937dff commit 5a5d290
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/data/fintype/basic.lean
Expand Up @@ -1515,7 +1515,7 @@ begin
intro; simp only [set.mem_to_finset, set.mem_compl_eq]; refl,
end

theorem card_subtype_mono (p q : α → Prop) (h : p ≤ q)
theorem fintype.card_subtype_mono (p q : α → Prop) (h : p ≤ q)
[fintype {x // p x}] [fintype {x // q x}] :
fintype.card {x // p x} ≤ fintype.card {x // q x} :=
fintype.card_le_of_embedding (subtype.imp_embedding _ _ h)
Expand Down

0 comments on commit 5a5d290

Please sign in to comment.