implication
Instances for implies
Implication →
is transitive. If P → Q
and Q → R
then P → R
.
not
false
eq
ne
and
or
xor
iff
iff P Q
, with notation P ↔ Q
, is the proposition asserting that P
and Q
are equivalent,
that is, have the same truth value.
Instances for iff
and simp rules
or simp rules
or resolution rulse
iff simp rules
implies simp rule
The existential quantifier.
To prove a goal of the form ⊢ ∃ x, p x
, you can provide a witness y
with the tactic existsi y
.
If you are working in a project that depends on mathlib, then we recommend the use
tactic
instead.
You'll then be left with the goal ⊢ p y
.
To extract a witness x
and proof hx : p x
from a hypothesis h : ∃ x, p x
,
use the tactic cases h with x hx
. See also the mathlib tactics obtain
and rcases
.
Instances for Exists
- exists_prop_decidable
- list.decidable_bex
- option.decidable_exists_mem
- bool.decidable_exists_bool
- nat.decidable_exists_lt
- nat.decidable_exists_le
- multiset.decidable_dexists_multiset
- finset.decidable_dexists_finset
- fintype.decidable_exists_fintype
- finset.decidable_exists_of_decidable_subsets
- finset.decidable_exists_of_decidable_ssubsets
- pnat.decidable_pred_exists_nat
exists unique
exists, forall, exists unique congruences
decidable
Equations
- decidable.to_bool p = h.cases_on (λ (h₁ : ¬p), bool.ff) (λ (h₂ : p), bool.tt)
Equations
Equations
Equations
- decidable.rec_on_true h₃ h₄ = h.rec_on (λ (h : ¬p), false.rec ((decidable.is_false h).rec_on h₂ h₁) _) (λ (h : p), h₄)
Equations
- decidable.rec_on_false h₃ h₄ = h.rec_on (λ (h : ¬p), h₄) (λ (h : p), false.rec ((decidable.is_true h).rec_on h₂ h₁) _)
Equations
- decidable_of_decidable_of_iff hp h = dite p (λ (hp : p), decidable.is_true _) (λ (hp : ¬p), decidable.is_false _)
Equations
Equations
- and.decidable = dite p (λ (hp : p), dite q (λ (hq : q), decidable.is_true _) (λ (hq : ¬q), decidable.is_false _)) (λ (hp : ¬p), decidable.is_false _)
Equations
- or.decidable = dite p (λ (hp : p), decidable.is_true _) (λ (hp : ¬p), dite q (λ (hq : q), decidable.is_true _) (λ (hq : ¬q), decidable.is_false _))
Equations
- not.decidable = dite p (λ (hp : p), decidable.is_false _) (λ (hp : ¬p), decidable.is_true hp)
Equations
- implies.decidable = dite p (λ (hp : p), dite q (λ (hq : q), decidable.is_true _) (λ (hq : ¬q), decidable.is_false _)) (λ (hp : ¬p), decidable.is_true _)
Equations
- iff.decidable = dite p (λ (hp : p), dite q (λ (hq : q), decidable.is_true _) (λ (hq : ¬q), decidable.is_false _)) (λ (hp : ¬p), dite q (λ (hq : q), decidable.is_false _) (λ (hq : ¬q), decidable.is_true _))
Equations
- xor.decidable = dite p (λ (hp : p), dite q (λ (hq : q), decidable.is_false _) (λ (hq : ¬q), decidable.is_true _)) (λ (hp : ¬p), dite q (λ (hq : q), decidable.is_true _) (λ (hq : ¬q), decidable.is_false _))
Equations
- exists_prop_decidable P = dite p (λ (h : p), decidable_of_decidable_of_iff (DP h) _) (λ (h : ¬p), decidable.is_false _)
Equations
- forall_prop_decidable P = dite p (λ (h : p), decidable_of_decidable_of_iff (DP h) _) (λ (h : ¬p), decidable.is_true _)
Equations
Equations
- decidable_eq_of_bool_pred h₁ h₂ = λ (x y : α), dite (p x y = bool.tt) (λ (hp : p x y = bool.tt), decidable.is_true _) (λ (hp : ¬p x y = bool.tt), decidable.is_false _)
inhabited
- default : α
Instances of this typeclass
- unique.inhabited
- prop.inhabited
- pi.inhabited
- bool.inhabited
- true.inhabited
- prod.inhabited
- nat.inhabited
- list.inhabited
- char.inhabited
- string.inhabited
- sum.inhabited_left
- sum.inhabited_right
- name.inhabited
- option.inhabited
- options.inhabited
- format.inhabited
- level.inhabited
- expr.inhabited
- environment.implicit_infer_kind.inhabited
- environment.inhabited
- local_context.inhabited
- occurrences.inhabited
- punit.inhabited
- json.inhabited
- sort.inhabited
- sort.inhabited'
- psum.inhabited_left
- psum.inhabited_right
- vm_decl_kind.inhabited
- vm_obj_kind.inhabited
- tactic.new_goals.inhabited
- tactic.transparency.inhabited
- tactic.apply_cfg.inhabited
- smt_pre_config.inhabited
- ematch_config.inhabited
- cc_config.inhabited
- smt_config.inhabited
- rsimp.config.inhabited
- tactic.dunfold_config.inhabited
- tactic.dsimp_config.inhabited
- tactic.unfold_proj_config.inhabited
- tactic.simp_intros_config.inhabited
- tactic.delta_config.inhabited
- tactic.simp_config.inhabited
- tactic.rewrite_cfg.inhabited
- interactive.loc.inhabited
- tactic.unfold_config.inhabited
- param_info.inhabited
- subsingleton_info.inhabited
- fun_info.inhabited
- format.color.inhabited
- pos.inhabited
- environment.projection_info.inhabited
- reducibility_hints.inhabited
- congr_arg_kind.inhabited
- ulift.inhabited
- plift.inhabited
- string_imp.inhabited
- string.iterator_imp.inhabited
- rbnode.color.inhabited
- ordering.inhabited
- unification_constraint.inhabited
- pprod.inhabited
- unification_hint.inhabited
- doc_category.inhabited
- tactic_doc_entry.inhabited
- bin_tree.inhabited
- unsigned.inhabited
- string.iterator.inhabited
- rbnode.inhabited
- rbtree.inhabited
- rbmap.inhabited
- binder_info.inhabited
- binder.inhabited
- tactic.goal.inhabited
- tactic.proof_state.inhabited
- to_additive.value_type.inhabited
- native.rb_set.inhabited
- native.rb_map.inhabited
- native.rb_lmap.inhabited
- name_set.inhabited
- name_map.inhabited
- lint_verbosity.inhabited
- tactic.rcases_patt.inhabited
- tactic.explode.status.inhabited
- tactic.explode.entries.inhabited
- auto.auto_config.inhabited
- auto.case_option.inhabited
- tactic.itauto.and_kind.inhabited
- tactic.itauto.prop.inhabited
- tactic.itauto.proof.inhabited
- norm_cast.label.inhabited
- norm_cast.norm_cast_cache.inhabited
- projection_data.inhabited
- simps_cfg.inhabited
- functor.const.inhabited
- functor.add_const.inhabited
- functor.comp.inhabited
- applicative_transformation.inhabited
- tactic.suggest.head_symbol_match.inhabited
- quot.inhabited
- quotient.inhabited
- trunc.inhabited
- fin.inhabited
- inhabited_fin_one_add
- units.inhabited
- add_units.inhabited
- equiv.inhabited'
- order_dual.inhabited
- as_linear_order.inhabited
- monoid.End.inhabited
- add_monoid.End.inhabited
- one_hom.inhabited
- zero_hom.inhabited
- mul_hom.inhabited
- add_hom.inhabited
- monoid_hom.inhabited
- add_monoid_hom.inhabited
- monoid_with_zero_hom.inhabited
- sigma.inhabited
- psigma.inhabited
- additive.inhabited
- multiplicative.inhabited
- mul_opposite.inhabited
- add_opposite.inhabited
- function.End.inhabited
- complementeds.inhabited
- with_bot.inhabited
- with_top.inhabited
- set.inhabited
- non_unital_ring_hom.inhabited
- ring_hom.inhabited
- mul_equiv.inhabited
- add_equiv.inhabited
- rel_embedding.inhabited
- rel_iso.inhabited
- tactic.interactive.mono_cfg.inhabited
- tactic.interactive.mono_selection.inhabited
- order_hom.inhabited
- with_one.inhabited
- with_zero.inhabited
- int.inhabited
- multiset.inhabited_multiset
- expr_lens.dir.inhabited
- tactic.interactive.rep_arity.inhabited
- finset.inhabited_finset
- pi.lex.inhabited
- pnat.inhabited
- rat.inhabited
- tactic.positivity.order_rel.inhabited
- top_hom.inhabited
- bot_hom.inhabited
- bounded_order_hom.inhabited
- sup_hom.inhabited
- inf_hom.inhabited
- sup_bot_hom.inhabited
- inf_top_hom.inhabited
- lattice_hom.inhabited
- bounded_lattice_hom.inhabited
- vector.inhabited
- sym.inhabited_sym
- sym.inhabited_sym'
- mul_aut.inhabited
- add_aut.inhabited
- tactic.abel.normalize_mode.inhabited
- ring_equiv.inhabited
- distrib_mul_action_hom.inhabited
- ring_aut.inhabited
- linear_map.inhabited
- associates.inhabited
- conj_classes.inhabited
- subsemigroup.inhabited
- add_subsemigroup.inhabited
- submonoid.inhabited
- add_submonoid.inhabited
- ulower.inhabited
- antisymmetrization.inhabited
- subgroup.inhabited
- add_subgroup.inhabited
- sub_mul_action.inhabited
- free_monoid.inhabited
- free_add_monoid.inhabited
- submodule.inhabited
- submodule.inhabited'
- set.finite.inhabited
- dfinsupp.inhabited
- finsupp.inhabited
- absolute_value.inhabited
- subsemiring.inhabited
- subring.inhabited
- alg_equiv.inhabited
- non_unital_alg_hom.inhabited
- tactic.tfae.arrow.inhabited
- part.inhabited
- omega_complete_partial_order.chain.inhabited
- omega_complete_partial_order.continuous_hom.inhabited
- monoid_algebra.inhabited
- add_monoid_algebra.inhabited
- polynomial.inhabited
- tactic.ring.normalize_mode.inhabited
- tactic.ring.ring_nf_cfg.inhabited
- linarith.ineq.inhabited
- linarith.comp.inhabited
- linarith.comp_source.inhabited
- prod.lex.inhabited
- pos_num.inhabited
- num.inhabited
- znum.inhabited
- tree.inhabited
- con.inhabited
- add_con.inhabited
- con.quotient.inhabited
- add_con.quotient.inhabited
- tensor_product.inhabited
- conj_act.inhabited
- Sup_hom.inhabited
- Inf_hom.inhabited
- frame_hom.inhabited
- complete_lattice_hom.inhabited
- set_semiring.inhabited
- enat.inhabited
- part_enat.inhabited
- cardinal.inhabited
- linear_pmap.inhabited
- quotient_group.has_quotient.quotient.inhabited
- quotient_add_group.has_quotient.quotient.inhabited
- submodule.quotient.has_quotient.quotient.inhabited
- basis.inhabited
- subalgebra.inhabited
- algebra.subalgebra.inhabited
- localization.inhabited
- add_localization.inhabited
- tactic.ring_exp.coeff.inhabited
- tactic.ring_exp.ex_type.inhabited
- zmod.inhabited
- restrict_scalars.inhabited
- unique_factorization_monoid.normalization_monoid.inhabited
- nat.primes.inhabited_primes
- cycle.inhabited
- mv_polynomial.inhabited
- ring_con.inhabited
- ring_con.quotient.inhabited
- ideal.quotient.inhabited
- local_ring.residue_field.inhabited
- direct_sum.inhabited
- self_adjoint.inhabited
- skew_adjoint.inhabited
- matrix.inhabited
- initial_seg.inhabited
- Well_order.inhabited
- ordinal.inhabited
- pequiv.inhabited
- composition_as_set.inhabited
- composition.inhabited
- nat.partition.inhabited
- multilinear_map.inhabited
- alternating_map.inhabited
- dmatrix.inhabited
- subfield.inhabited
- intermediate_field.alg_hom.inhabited
- perfect_closure.inhabited
- free_algebra.pre.inhabited
- free_algebra.inhabited
- adjoin_root.inhabited
- intermediate_field.inhabited
- intermediate_field.lifts.inhabited
- abelianization.inhabited
- polynomial.splitting_field_aux.inhabited
- polynomial.splitting_field.inhabited
- lift.subfield_with_hom.inhabited
- galois_field.inhabited
- filter.inhabited_mem
- filter.inhabited
- filter_basis.inhabited
- filter.nat.inhabited_countable_filter_basis
- tactic.decl_reducibility.inhabited
- ultrafilter.inhabited
- inhabited_topological_space
- cofinite_topology.inhabited
- upper_set.inhabited
- lower_set.inhabited
- compact_exhaustion.inhabited
- connected_components.inhabited
- separation_quotient.inhabited
- inhabited_uniform_space
- inhabited_uniform_space_core
- uniform_space.separation_quotient.inhabited
- continuous_map.inhabited
- group_topology.inhabited
- add_group_topology.inhabited
- ring_topology.inhabited
- nonneg.inhabited
- cau_seq.inhabited
- cau_seq.completion.Cauchy.inhabited
- real.inhabited
- nnreal.inhabited
- ennreal.inhabited
- Cauchy.inhabited
- uniform_space.completion.inhabited
- uniform_space.completion.abstract_completion.inhabited
- complex.inhabited
- group_seminorm.inhabited
- add_group_seminorm.inhabited
- nonarch_add_group_seminorm.inhabited
- add_group_norm.inhabited
- group_norm.inhabited
- nonarch_add_group_norm.inhabited
- locally_bounded_map.inhabited
- normed_add_group_hom.inhabited
- continuous_linear_map.inhabited
- linear_isometry.inhabited
- linear_isometry_equiv.inhabited
- unitary.inhabited
- non_unital_star_alg_hom.inhabited
- star_alg_hom.inhabited
- star_alg_equiv.inhabited
- star_subalgebra.inhabited
- list.tprod.inhabited
- measurable_space.inhabited
- measurable_space.dynkin_system.inhabited
- measure_theory.outer_measure.inhabited
- measurable_equiv.inhabited
- measure_theory.null_measurable_space.inhabited
- measure_theory.measure.inhabited
- derive_fintype.finset_above.inhabited
- sign_type.inhabited
- ereal.inhabited
- measure_theory.simple_func.inhabited
- cocompact_map.inhabited
- stieltjes_function.inhabited
- topological_space.opens.inhabited
- topological_space.open_nhds_of.inhabited
- topological_space.closeds.inhabited
- topological_space.clopens.inhabited
- topological_space.compacts.inhabited
- topological_space.nonempty_compacts.inhabited
- topological_space.positive_compacts.inhabited
- topological_space.compact_opens.inhabited
- measure_theory.content.inhabited
- affine_map.inhabited
- affine_subspace.inhabited
- module.dual.inhabited
- bilin_form.inhabited
- closure_operator.inhabited
- lower_adjoint.inhabited
- affine.simplex.inhabited
- affine_basis.inhabited
- zeroth_homotopy.inhabited
- affine_isometry.inhabited
- affine_isometry_equiv.inhabited
- local_equiv.inhabited
- local_equiv.inhabited_of_empty
- seminorm.inhabited
- group_filter_basis.inhabited
- add_group_filter_basis.inhabited
- module_filter_basis.inhabited
- continuous_multilinear_map.inhabited
- continuous_linear_map.nonlinear_right_inverse.inhabited
- composition_series.inhabited
- add_circle.inhabited
- real.angle.inhabited
- pi_Lp.inhabited
- orthonormal_basis.inhabited
- box_integral.box.inhabited
- box_integral.prepartition.inhabited
- box_integral.tagged_prepartition.inhabited
- box_integral.integration_params.inhabited
- box_integral.box_additive_map.inhabited
- filter.product.inhabited
- filter.germ.inhabited
- urysohns.CU.inhabited
- bounded_continuous_function.inhabited
- measure_theory.ae_eq_fun.inhabited
- formal_multilinear_series.inhabited
- matrix.special_linear_group.inhabited
- convex_cone.inhabited
- weak_dual.inhabited
- normed_space.dual.inhabited
- mv_power_series.inhabited
- power_series.inhabited
- hahn_series.inhabited
- hahn_series.summable_family.inhabited
- ratfunc.inhabited
- open_subgroup.inhabited
- open_add_subgroup.inhabited
- free_group.inhabited
- free_add_group.inhabited
- free_abelian_group.inhabited
- free_ring.inhabited
- free_comm_ring.inhabited
- module.direct_limit.inhabited
- add_comm_group.direct_limit.inhabited
- ring.direct_limit.inhabited
- algebraic_closure.adjoin_monic.inhabited
- algebraic_closure.step.inhabited
- algebraic_closure.inhabited
- mv_polynomial.R.inhabited
- opposite.inhabited
- prefunctor.inhabited
- lazy_list.inhabited
- slim_check.no_shrink.inhabited
- slim_check.small.inhabited
- slim_check.large.inhabited
- slim_check.test_result.inhabited
- slim_check.slim_check_cfg.inhabited
- slim_check.use_has_to_string.inhabited
- d_array.inhabited
- array.inhabited
- buffer.inhabited
- parser.inhabited
- polyrith.poly.inhabited
- polyrith.sage_json_success.inhabited
- polyrith.sage_json_failure.inhabited
- tactic.eliminate.generalization_mode.inhabited
- nzsnum.inhabited
- snum.inhabited
- tactic.ring2.csring_expr.inhabited
- tactic.ring2.horner_expr.inhabited
- omega.term.inhabited
- omega.ee.inhabited
- omega.ee_state.inhabited
- omega.int.preterm.inhabited
- omega.int.preform.inhabited
- omega.nat.preterm.inhabited
- omega.nat.preform.inhabited
- category_theory.functor.inhabited
- category_theory.nat_trans.inhabited
- category_theory.iso.inhabited
- category_theory.equivalence.inhabited
- quiver.wide_subquiver.inhabited
- quiver.labelling.inhabited
- quiver.path.inhabited
- quiver.weakly_connected_component.inhabited
- category_theory.comma.inhabited
- category_theory.comma_morphism.inhabited
- category_theory.arrow.inhabited
- category_theory.adjunction.inhabited
- category_theory.discrete.inhabited
- category_theory.limits.inhabited_cone
- category_theory.limits.inhabited_cocone
- category_theory.limits.inhabited_cone_morphism
- category_theory.limits.inhabited_cocone_morphism
- category_theory.ulift_hom.inhabited
- category_theory.as_small.inhabited
- category_theory.limits.wide_pullback_shape.inhabited
- category_theory.limits.wide_pushout_shape.inhabited
- category_theory.limits.wide_pullback_shape.hom.inhabited
- category_theory.limits.wide_pushout_shape.hom.inhabited
- category_theory.Cat.inhabited
- category_theory.skeleton.inhabited
- category_theory.inhabited_thin_skeleton
- category_theory.thin_skeleton.is_skeleton_of_inhabited
- category_theory.over.inhabited
- category_theory.under.inhabited
- category_theory.limits.walking_pair.inhabited
- tactic.rewrite_search.side.inhabited
- tactic.rewrite_search.dir_pair.inhabited
- tactic.rewrite_search.using_conv.splice_result.inhabited
- side.inhabited
- measure_theory.vector_measure.inhabited
- measure_theory.jordan_decomposition.inhabited
- measure_theory.filtration.inhabited
- metric.inhabited_left
- metric.inhabited_right
- metric.inductive_limit.inhabited
- pmf.inhabited
- representation.as_module.inhabited
- Mon.inhabited
- AddMon.inhabited
- CommMon.inhabited
- AddCommMon.inhabited
- category_theory.End.inhabited
- category_theory.Aut.inhabited
- Group.inhabited
- AddGroup.inhabited
- CommGroup.inhabited
- AddCommGroup.inhabited
- quiver.single_obj.inhabited
- category_theory.inhabited_liftable_cone
- category_theory.inhabited_liftable_cocone
- category_theory.inhabited_lifts_to_limit
- category_theory.inhabited_lifts_to_colimit
- category_theory.lax_monoidal_functor.inhabited
- category_theory.monoidal_functor.inhabited
- category_theory.free_monoidal_category.inhabited
- hom_rel.inhabited
- category_theory.quotient.inhabited
- category_theory.quotient.hom.inhabited
- category_theory.paths.inhabited
- category_theory.prelax_functor.inhabited
- category_theory.oplax_functor.inhabited
- category_theory.pseudofunctor.inhabited
- category_theory.free_bicategory.inhabited
- category_theory.free_bicategory.hom.inhabited
- category_theory.locally_discrete.inhabited
- category_theory.monoidal_nat_trans.inhabited
- category_theory.lax_braided_functor.inhabited
- category_theory.braided_functor.inhabited
- category_theory.monoidal.transported.inhabited
- category_theory.limits.walking_parallel_pair.inhabited
- category_theory.limits.walking_parallel_pair_hom.inhabited
- category_theory.limits.mono_factorisation.inhabited
- category_theory.limits.is_image.inhabited
- category_theory.limits.image_factorisation.inhabited
- category_theory.limits.inhabited_image_map
- category_theory.limits.strong_epi_mono_factorisation_inhabited
- category_theory.limits.types.image.inhabited
- category_theory.is_split_coequalizer.inhabited
- Action.inhabited'
- Action.inhabited
- Action.hom.inhabited
- Module.inhabited
- category_theory.mono_over.inhabited
- category_theory.subobject.inhabited
- Module.colimits.prequotient.inhabited
- Module.colimits.colimit_type.inhabited
- fgModule.inhabited
- category_theory.inhabited_graded_object
- homological_complex.hom.inhabited
- homological_complex.inhabited
- Fintype.inhabited
- Fintype.skeleton.inhabited
- Preord.inhabited
- PartOrd.inhabited
- FinPartOrd.inhabited
- Lat.inhabited
- LinOrd.inhabited
- NonemptyFinLinOrd.inhabited
- simplex_category.inhabited
- simplex_category.truncated.inhabited
- category_theory.idempotents.karoubi.hom.inhabited
- Top.inhabited
- category_theory.limits.walking_multicospan.inhabited
- category_theory.limits.walking_multicospan.hom.inhabited
- category_theory.limits.walking_multispan.inhabited
- category_theory.limits.walking_multispan.hom.inhabited
- sSet.inhabited
- sSet.truncated.inhabited
- homotopy_equiv.inhabited
- homotopy_category.inhabited
- category_theory.abelian.pseudoelement.inhabited
- besicovitch.satellite_config.inhabited
- besicovitch.ball_package.inhabited
- besicovitch.tau_package.inhabited
- measure_theory.finite_measure.inhabited
- measure_theory.probability_measure.inhabited
- category_theory.monad_hom.inhabited
- category_theory.comonad_hom.inhabited
- category_theory.monad.inhabited
- category_theory.comonad.inhabited
- category_theory.monad.algebra.hom.inhabited
- category_theory.monad.algebra.inhabited
- Meas.inhabited
- continuous_affine_map.inhabited
- stone_cech.inhabited
- alexandroff.inhabited
- bump_covering.inhabited
- partition_of_unity.inhabited
- rel.inhabited
- pfun.inhabited
- bundle.total_space.inhabited
- locally_constant.inhabited
- discrete_quotient.inhabited
- discrete_quotient.inhabited_quotient
- triv_sq_zero_ext.inhabited
- spectral_map.inhabited
- clopen_upper_set.inhabited
- Gromov_Hausdorff.GH_space.inhabited
- Gromov_Hausdorff.aux_gluing_struct.inhabited
- dilation.inhabited
- vector_bundle_core.inhabited
- continuous_map.homotopy.inhabited
- continuous_map.homotopy_with.inhabited
- path.homotopic.quotient.inhabited
- category_theory.Groupoid.inhabited
- fundamental_groupoid.inhabited
- fundamental_group.inhabited
- loop_space.inhabited
- gen_loop.inhabited
- homotopy_group.inhabited
- continuous_map.homotopy_equiv.inhabited
- with_lower_topology.inhabited
- continuous_order_hom.inhabited
- pseudo_epimorphism.inhabited
- esakia_hom.inhabited
- continuous_open_map.inhabited
- compare_reals.Q.inhabited
- compare_reals.Bourbakiℝ.inhabited
- UniformSpace.inhabited
- CpltSepUniformSpace.inhabited
- SemiRing.inhabited
- Ring.inhabited
- CommSemiRing.inhabited
- CommRing.inhabited
- TopCommRing.inhabited
- Born.inhabited
- CompHaus.inhabited
- Frm.inhabited
- Locale.inhabited
- category_theory.kleisli.inhabited
- category_theory.cokleisli.inhabited
- category_theory.Kleisli.inhabited
- category_theory.Kleisli.mk.inhabited
- Profinite.inhabited
- Compactum.inhabited
- topological_space.open_nhds.inhabited
- continuous_monoid_hom.inhabited
- continuous_add_monoid_hom.inhabited
- pontryagin_dual.inhabited
- derivation.inhabited
- zero_at_infty_continuous_map.inhabited
- category_theory.presieve.inhabited
- category_theory.sieve.sieve_inhabited
- category_theory.grothendieck_topology.inhabited
- category_theory.grothendieck_topology.cover.inhabited
- category_theory.pretopology.inhabited
- category_theory.presieve.family_of_elements.inhabited
- category_theory.equalizer.first_obj.inhabited
- category_theory.equalizer.sieve.second_obj.inhabited
- category_theory.equalizer.presieve.second_obj.inhabited
- category_theory.SheafOfTypes.hom.inhabited
- category_theory.SheafOfTypes.inhabited
- category_theory.Sheaf.hom.inhabited
- category_theory.Sheaf.inhabited
- Top.sheaf_inhabited
- category_theory.bicone.inhabited
- category_theory.bicone_hom.inhabited
- Top.presheaf.sheaf_condition.opens_le_cover.inhabited
- category_theory.pairwise.pairwise_inhabited
- category_theory.pairwise.hom_inhabited
- CommRing.colimits.prequotient.inhabited
- CommRing.colimits.colimit_type.inhabited
- Top.presheaf.submonoid_presheaf.inhabited
- Top.inhabited_prelocal_predicate
- Top.inhabited_local_predicate
- category_theory.subterminals.inhabited
- category_theory.grothendieck.hom.inhabited
- category_theory.with_terminal.inhabited
- category_theory.with_initial.inhabited
- category_theory.is_kernel_pair.inhabited
- category_theory.morphism_property.inhabited
- semidirect_product.inhabited
- category_theory.action_category.inhabited
- category_theory.sigma.sigma_hom.inhabited
- category_theory.connected_components.inhabited
- category_theory.component.inhabited
- category_theory.oplax_nat_trans.inhabited
- category_theory.oplax_nat_trans.modification.inhabited
- category_theory.End_monoidal.inhabited
- category_theory.monoidal_single_obj.inhabited
- category_theory.endofunctor.algebra.inhabited
- category_theory.endofunctor.algebra.hom.inhabited
- category_theory.endofunctor.coalgebra.inhabited
- category_theory.endofunctor.coalgebra.hom.inhabited
- category_theory.subgroupoid.inhabited
- category_theory.limits.diagram_of_cones_inhabited
- category_theory.parallel_pair_inhabited
- category_theory.limits.walking_parallel_family.inhabited
- category_theory.limits.walking_parallel_family.hom.inhabited
- category_theory.Mat_.quiver.hom.inhabited
- category_theory.Mat_.inhabited
- category_theory.Mat.inhabited
- category_theory.Mat.quiver.hom.inhabited
- Pointed.inhabited
- Pointed.hom.inhabited
- Bipointed.inhabited
- Bipointed.hom.inhabited
- two_pointing.inhabited
- Twop.inhabited
- category_theory.Quiv.inhabited
- category_theory.Rel.inhabited
- PartialFun.inhabited
- category_theory.localization.strict_universal_property_fixed_target.inhabited
- category_theory.pretriangulated.triangle.inhabited
- category_theory.pretriangulated.triangle_morphism.inhabited
- Mon_.inhabited
- Mon_.hom_inhabited
- Bimod.hom_inhabited
- Bimod.inhabited
- Mod_.hom_inhabited
- Mod_.inhabited
- CommMon_.inhabited
- Mon_Type_inhabited
- CommMon_Type_inhabited
- Algebra.inhabited
- category_theory.enriched_functor.inhabited
- flow.inhabited
- circle_deg1_lift.inhabited
- stream.inhabited
- fin2.inhabited
- typevec.inhabited
- typevec.arrow.inhabited
- typevec.last.inhabited
- typevec.curry.inhabited
- schwartz_map.inhabited
- cont_diff_bump.inhabited
- quaternion_algebra.inhabited
- quaternion.inhabited
- hilbert_basis.inhabited
- polynomial_module.inhabited
- picard_lindelof.inhabited
- picard_lindelof.fun_space.inhabited
- enorm.inhabited
- double_centralizer.inhabited
- ring_seminorm.inhabited
- ring_norm.inhabited
- mul_ring_seminorm.inhabited
- mul_ring_norm.inhabited
- SemiNormedGroup.inhabited
- SemiNormedGroup₁.inhabited
- upper_half_plane.inhabited
- structure_groupoid.inhabited
- pregroupoid.inhabited
- model_prod_inhabited
- model_pi_inhabited
- tangent_space.inhabited
- cont_mdiff_map.inhabited
- complex.unit_disc.inhabited
- convex_body.inhabited
- geometry.simplicial_complex.inhabited
- proper_cone.inhabited
- ideal.cotangent.inhabited
- perfection.ring.perfection.inhabited
- ring_invo.inhabited
- fractional_ideal.inhabited
- class_group.inhabited
- ideal.filtration.inhabited
- non_unital_subsemiring.inhabited
- graded_monoid.inhabited
- homogeneous_ideal.inhabited
- ore_localization.inhabited
- witt_vector.inhabited
- witt_vector.is_poly.inhabited
- witt_vector.is_poly₂.inhabited
- truncated_witt_vector.inhabited
- padic.inhabited
- padic_int.inhabited
- valuation_ring.value_group.inhabited
- valuation_subring.inhabited
- valuation_subring.inhabited_value_group
- is_dedekind_domain.height_one_spectrum.adic_completion.inhabited
- is_dedekind_domain.height_one_spectrum.adic_completion_integers.inhabited
- dedekind_domain.finite_integral_adeles.inhabited
- dedekind_domain.prod_adic_completions.inhabited
- lie_hom.inhabited
- lie_equiv.inhabited
- lie_module_hom.inhabited
- lie_module_equiv.inhabited
- lie_subalgebra.inhabited
- lie_submodule.inhabited
- nat.arithmetic_function.inhabited
- nonempty_interval.inhabited
- interval.inhabited
- order.ideal.inhabited
- order.cofinal.inhabited
- order.pfilter.inhabited
- concept.inhabited
- order.partial_iso.inhabited
- well_order_extension.inhabited
- linear_extension.inhabited
- finpartition.inhabited
- heyting_hom.inhabited
- coheyting_hom.inhabited
- biheyting_hom.inhabited
- heyting.regular.inhabited
- BddOrd.inhabited
- SemilatSup.inhabited
- SemilatInf.inhabited
- BddLat.inhabited
- DistLat.inhabited
- BddDistLat.inhabited
- HeytAlg.inhabited
- BoolAlg.inhabited
- FinBddDistLat.inhabited
- FinBoolAlg.inhabited
- CompleteLat.inhabited
- ωCPO.inhabited
- simplicial_object.splitting.index_set.inhabited
- computation.inhabited
- stream.seq.inhabited
- stream.seq1.inhabited
- generalized_continued_fraction.pair.inhabited
- generalized_continued_fraction.inhabited
- simple_continued_fraction.inhabited
- continued_fraction.inhabited
- generalized_continued_fraction.int_fract_pair.inhabited
- zsqrtd.inhabited
- pell.solution₁.inhabited
- mul_char.inhabited
- cyclotomic_field.inhabited
- cyclotomic_ring.inhabited
- add_char.inhabited
- lucas_lehmer.X.inhabited
- function_field.Fqt_infty.inhabited
- vector3.inhabited
- poly.inhabited
- slash_invariant_form.inhabited
- modular_form.inhabited
- cusp_form.inhabited
- absolute_value.is_admissible.inhabited
- smooth_bump_function.inhabited
- smooth_monoid_morphism.inhabited
- smooth_add_monoid_morphism.inhabited
- smooth_partition_of_unity.inhabited
- euclidean_half_space.inhabited
- euclidean_quadrant.inhabited
- pointed_smooth_map.inhabited
- cont_mdiff_section.inhabited
- left_invariant_derivation.inhabited
- affine.simplex.points_with_circumcenter_index_inhabited
- lists'.inhabited
- lists.inhabited
- finsets.inhabited
- pgame.inhabited
- pgame.relabelling.inhabited
- game.inhabited
- pgame.inv_ty.inhabited
- nat_ordinal.inhabited
- order_monoid_hom.inhabited
- order_add_monoid_hom.inhabited
- order_monoid_with_zero_hom.inhabited
- surreal.inhabited
- arity.arity.inhabited
- pSet.inhabited
- pSet.type.inhabited
- pSet.resp.inhabited
- Set.inhabited
- Class.inhabited
- onote.inhabited
- nonote.inhabited
- pgame.domineering.board.inhabited
- ring_quot.inhabited
- shelf_hom.inhabited
- rack.pre_envel_group.inhabited
- rack.pre_envel_group_rel'.inhabited
- rack.envel_group.inhabited
- free_magma.inhabited
- free_add_magma.inhabited
- magma.assoc_quotient.inhabited
- add_magma.free_add_semigroup.inhabited
- free_semigroup.inhabited
- free_add_semigroup.inhabited
- cubic.inhabited
- linear_recurrence.inhabited
- quaternion_algebra.basis.inhabited
- sym_alg.inhabited
- as_boolalg.inhabited
- as_boolring.inhabited
- tropical.inhabited
- module.Baer.extension_of.inhabited
- local_cohomology.self_le_radical.inhabited
- lie_submodule.quotient.inhabited
- lie_algebra.commutator_ring.inhabited
- tensor_algebra.inhabited
- universal_enveloping_algebra.inhabited
- free_lie_algebra.inhabited
- cartan_matrix.generators.inhabited
- matrix.to_lie_algebra.inhabited
- order_ring_hom.inhabited
- order_ring_iso.inhabited
- freiman_hom.inhabited
- add_freiman_hom.inhabited
- centroid_hom.inhabited
- GroupWithZero.inhabited
- BoolRing.inhabited
- AddCommGroup.colimits.prequotient.inhabited
- AddCommGroup.colimits.colimit_type.inhabited
- Mon.colimits.prequotient.inhabited
- Mon.colimits.colimit_type.inhabited
- Magma.inhabited
- AddMagma.inhabited
- Semigroup.inhabited
- AddSemigroup.inhabited
- unitization.inhabited
- pi_tensor_product.inhabited
- quadratic_form.inhabited
- clifford_algebra.inhabited
- clifford_algebra.even_hom.inhabited
- module.End.eigenvalues.inhabited
- projectivization.subspace.subspace_inhabited
- language.inhabited
- DFA.inhabited
- NFA.inhabited
- ε_NFA.inhabited
- regular_expression.inhabited
- nat.partrec.code.inhabited
- turing.list_blank.inhabited
- turing.pointed_map.inhabited
- turing.tape.inhabited
- turing.dir.inhabited
- turing.TM0.stmt.inhabited
- turing.TM0.machine.inhabited
- turing.TM0.cfg.inhabited
- turing.TM1.stmt.inhabited
- turing.TM1.cfg.inhabited
- turing.TM1to0.Λ'.inhabited
- turing.TM1to1.Λ'.inhabited
- turing.TM0to1.Λ'.inhabited
- turing.TM2.stmt.inhabited
- turing.TM2.cfg.inhabited
- turing.TM2to1.Γ'.inhabited
- turing.TM2to1.st_act.inhabited
- turing.TM2to1.Λ'.inhabited
- turing.to_partrec.code.inhabited
- turing.to_partrec.cont.inhabited
- turing.to_partrec.cfg.inhabited
- turing.partrec_to_TM2.Γ'.inhabited
- turing.partrec_to_TM2.K'.inhabited
- turing.partrec_to_TM2.cont'.inhabited
- turing.partrec_to_TM2.Λ'.inhabited
- turing.partrec_to_TM2.stmt'.inhabited
- turing.partrec_to_TM2.cfg'.inhabited
- computability.inhabited_Γ'
- computability.inhabited_fin_encoding
- computability.inhabited_encoding
- turing.fin_tm2.σ.inhabited
- turing.fin_tm2.stmt.inhabited
- turing.fin_tm2.inhabited_cfg
- turing.inhabited_fin_tm2
- turing.inhabited_tm2_computable_in_poly_time
- turing.inhabited_tm2_outputs_in_time
- turing.inhabited_tm2_outputs
- turing.inhabited_evals_to_in_time
- turing.inhabited_tm2_evals_to
- turing.inhabited_tm2_computable_in_time
- turing.inhabited_tm2_computable
- turing.inhabited_tm2_computable_aux
- many_one_degree.inhabited
- slim_check.total_function.inhabited
- slim_check.injective_function.inhabited
- combinatorics.line.inhabited
- combinatorics.line.almost_mono.inhabited
- combinatorics.line.color_focused.inhabited
- finset.colex.inhabited
- configuration.dual.inhabited
- nnrat.inhabited
- simple_graph.inhabited
- indexed_partition.inhabited
- indexed_partition.quotient.inhabited
- simple_graph.partition.inhabited
- simple_graph.subgraph.subgraph_inhabited
- simple_graph.walk.inhabited
- simple_graph.connected_component.inhabited
- young_diagram.inhabited
- ssyt.inhabited
- semiquot.inhabited
- erased.inhabited
- bucket_array.inhabited
- hash_map.inhabited
- alist.inhabited
- finmap.inhabited
- holor.inhabited
- W_type.inhabited
- W_type.nat_α.inhabited
- W_type.nat_β.inhabited
- W_type.list_α.inhabited
- W_type.list_β.inhabited
- pfunctor.inhabited
- pfunctor.obj.inhabited
- pfunctor.Idx.inhabited
- mvpfunctor.inhabited
- mvpfunctor.obj.inhabited
- pfunctor.approx.cofix_a.inhabited
- pfunctor.approx.path.inhabited
- pfunctor.M.inhabited
- pfunctor.M_intl.inhabited
- mvpfunctor.M.path.inhabited
- mvpfunctor.inhabited_M
- mvqpf.cofix.inhabited
- mvqpf.prj.inhabited
- mvqpf.comp.inhabited
- mvqpf.quot1.inhabited
- mvpfunctor.W_path.inhabited
- mvqpf.const.inhabited
- mvqpf.sigma.inhabited
- mvqpf.pi.inhabited
- qpf.cofix.inhabited
- stream.wseq.inhabited
- hyperreal.inhabited
- cfilter.inhabited
- filter.realizer.realizer.inhabited
- ctop.inhabited
- ctop.realizer.inhabited
- compact.realizer.inhabited
- prime_multiset.inhabited
- pnat.xgcd_type.inhabited
- ordnode.inhabited
- ordset.inhabited
- dlist.inhabited
- fp.rmode.inhabited
- fp.float.inhabited
- hamming.inhabited
- first_order.sequence₂.inhabited₀
- first_order.sequence₂.inhabited₁
- first_order.sequence₂.inhabited₂
- first_order.language.inhabited
- first_order.language.hom.inhabited
- first_order.language.embedding.inhabited
- first_order.language.equiv.inhabited
- first_order.language.Lhom.inhabited
- first_order.language.Lequiv.inhabited
- first_order.language.term.inhabited_of_var
- first_order.language.term.inhabited_of_constant
- first_order.language.bounded_formula.inhabited
- first_order.language.substructure.inhabited
- first_order.language.direct_limit.inhabited
- first_order.language.elementary_embedding.inhabited
- first_order.language.elementary_substructure.inhabited
- first_order.language.Theory.Model.inhabited
- first_order.language.definable_set.inhabited
- algebraic_geometry.PresheafedSpace.inhabited
- algebraic_geometry.PresheafedSpace.hom_inhabited
- algebraic_geometry.SheafedSpace.inhabited
- algebraic_geometry.LocallyRingedSpace.hom.inhabited
- algebraic_geometry.structure_sheaf.localizations.inhabited
- algebraic_geometry.Scheme.inhabited
- algebraic_geometry.Scheme.open_cover.inhabited
- weierstrass_curve.inhabited
- weierstrass_curve.coordinate_ring.inhabited
- elliptic_curve.inhabited
- weierstrass_curve.point.inhabited
- algebraic_geometry.affine_target_morphism_property.inhabited
- sylow.inhabited
- subgroup.left_transversals.inhabited
- add_subgroup.left_transversals.inhabited
- subgroup.right_transversals.inhabited
- add_subgroup.right_transversals.inhabited
- free_product.inhabited
- free_product.word.inhabited
- free_product.word.pair.inhabited
- subgroup.quotient_diff.inhabited
- presented_group.inhabited
- doset.quotient.inhabited
- dihedral_group.inhabited
- quaternion_group.inhabited
- counterexample.int_with_epsilon.inhabited
- counterexample.F.inhabited
- counterexample.from_Bhavik.inhabited_K
- counterexample.ex_L.inhabited
- counterexample.foo.inhabited
- counterexample.discrete_copy.inhabited
- counterexample.phillips_1940.bounded_additive_measure.inhabited
- arithcc.expr.inhabited
- arithcc.instruction.inhabited
- arithcc.state.inhabited
- sensitivity.Q.inhabited
- miu.miu_atom_inhabited
Instances of other typeclasses for inhabited
- inhabited.has_sizeof_inst
Equations
- prop.inhabited = {default := true}
Equations
- pi.inhabited α = {default := λ (a : α), inhabited.default}
Equations
Equations
Instances of this typeclass
- has_zero.nonempty
- has_one.nonempty
- has_Inf_to_nonempty
- has_Sup_to_nonempty
- irreducible_space.to_nonempty
- connected_space.to_nonempty
- has_top_nonempty
- has_bot_nonempty
- add_torsor.nonempty
- category_theory.is_connected.is_nonempty
- nontrivial.to_nonempty
- nonempty_of_inhabited
- prod.nonempty
- pi.nonempty
- order_dual.nonempty
- nonempty_lt
- nonempty_gt
- set.univ.nonempty
- set.has_insert.insert.nonempty
- set.image.nonempty
- set.range.nonempty
- set.nonempty_Ici_subtype
- set.nonempty_Iic_subtype
- set.nonempty_Ioi_subtype
- set.nonempty_Iio_subtype
- plift.nonempty
- ulift.nonempty
- finset.has_insert.insert.nonempty
- nonempty_equiv_of_countable
- commutator_set.nonempty
- module.free.choose_basis_index.nonempty
- is_well_order.subtype_nonempty
- cardinal.nonempty_out_aleph
- filter_basis.nonempty_sets
- ultrafilter.nonempty
- separation_quotient.nonempty
- uniform_fun.nonempty
- uniform_on_fun.nonempty
- Cauchy.nonempty
- matrix.transvection_struct.nonempty
- topological_space.nonempty_compacts.to_nonempty
- topological_space.positive_compacts.nonempty'
- affine_map.nonempty
- ray_vector.nonempty
- module.ray.nonempty
- affine_span.nonempty
- affine.simplex.nonempty
- unit_interval.nonempty
- quiver.push.nonempty
- nonempty_fin_lin_ord.nonempty
- sSet.augmented.standard_simplex.nonempty_extra_degeneracy_standard_simplex
- bundle.pullback.nonempty
- discrete_quotient.nonempty
- Gromov_Hausdorff.rep_GH_space_nonempty
- with_lower_topology.nonempty
- category_theory.nonempty_hom_of_connected_groupoid
- category_theory.functor.final.category_theory.structured_arrow.nonempty
- category_theory.functor.initial.category_theory.costructured_arrow.nonempty
- Top.presheaf.sheaf_condition.category_theory.structured_arrow.nonempty
- category_theory.grothendieck_topology.subpresheaf.nonempty
- category_theory.action_category.nonempty
- category_theory.component.nonempty
- category_theory.groupoid.free.category_theory.free_groupoid.nonempty
- two_pointing.nonempty
- category_theory.triangulated.octahedron.nonempty
- weak_dual.character_space.nonempty
- abs_convex_open_sets.nonempty
- kaehler_differential.nonempty
- prime_spectrum.nonempty
- maximal_spectrum.nonempty
- nonempty_interval.nonempty
- set.subchain.nonempty
- number_field.embeddings.ring_hom.nonempty
- number_field.infinite_place.nonempty
- euclidean_geometry.sphere.nonempty
- lie_algebra.commutator_ring.nonempty
- projectivization.nonempty
- quiver.rooted_connected.nonempty_path
- simple_graph.nonempty_dart_top
- simple_graph.nonempty_singleton_subgraph_verts
- simple_graph.nonempty_subgraph_of_adj_verts
- locally_finite.realizer.nonempty
- first_order.language.elementary_substructure.nonempty
- first_order.language.Theory.Model.nonempty'
- first_order.language.Theory.Model.nonempty
- first_order.language.ultraproduct.product.nonempty
- first_order.language.Theory.complete_type.nonempty
- algebraic_geometry.is_integral.nonempty
- sylow.nonempty
subsingleton
Instances of this typeclass
- is_empty.subsingleton
- unique.subsingleton
- char_p.subsingleton
- category_theory.quiver.is_thin
- subsingleton_prop
- decidable.subsingleton
- pi.subsingleton
- punit.subsingleton
- empty.subsingleton
- subsingleton.prod
- subtype.subsingleton
- subsingleton_pempty
- quot.subsingleton
- quotient.subsingleton
- trunc.subsingleton
- unique.subsingleton_unique
- equiv.equiv_subsingleton_cod
- equiv.equiv_subsingleton_dom
- order_dual.subsingleton
- mul_opposite.subsingleton
- add_opposite.subsingleton
- invertible.subsingleton
- set.subsingleton_coe_of_subsingleton
- ring_hom.int.subsingleton_ring_hom
- fin.order_iso_subsingleton
- fin.order_iso_subsingleton'
- plift.subsingleton
- ulift.subsingleton
- fintype.subsingleton
- rat.subsingleton_ring_hom
- vector.zero_subsingleton
- sym.subsingleton
- subsingleton_rat_module
- subsingleton_gcd_monoid_of_unique_units
- subsingleton_normalized_gcd_monoid_of_unique_units
- subsingleton_fin_zero
- subsingleton_fin_one
- nat_algebra_subsingleton
- algebra_rat_subsingleton
- int_algebra_subsingleton
- locally_finite_order.subsingleton
- locally_finite_order_top.subsingleton
- locally_finite_order_bot.subsingleton
- order.succ_order.subsingleton
- order.pred_order.subsingleton
- subalgebra.subsingleton_of_subsingleton
- alg_hom.subsingleton
- alg_equiv.subsingleton_left
- alg_equiv.subsingleton_right
- matrix.subsingleton
- matrix.subsingleton_of_empty_left
- matrix.subsingleton_of_empty_right
- initial_seg.subsingleton_of_trichotomous_of_irrefl
- initial_seg.subsingleton
- principal_seg.subsingleton
- dmatrix.subsingleton
- dmatrix.subsingleton_of_empty_left
- dmatrix.subsingleton_of_empty_right
- zmod.subsingleton_units
- zmod.subsingleton_ring_hom
- zmod.subsingleton_ring_equiv
- zmod.algebra.subsingleton
- separation_quotient.subsingleton
- measure_theory.null_measurable_space.subsingleton
- measure_theory.measure.subsingleton
- direct_sum.decomposition.subsingleton
- continuous_map.subsingleton_subalgebra
- hahn_series.subsingleton
- ratfunc.subsingleton
- category_theory.subsingleton_of_unop
- category_theory.comm_sq.subsingleton_lift_struct_of_epi
- category_theory.comm_sq.subsingleton_lift_struct_of_mono
- category_theory.discrete.subsingleton
- category_theory.limits.is_limit.subsingleton
- category_theory.limits.is_colimit.subsingleton
- category_theory.functor_thin
- category_theory.subsingleton_iso
- category_theory.limits.wide_pullback_shape.subsingleton_hom
- category_theory.limits.wide_pushout_shape.subsingleton_hom
- category_theory.thin_skeleton.thin
- category_theory.limits.walking_cospan.quiver.hom.subsingleton
- category_theory.limits.walking_span.quiver.hom.subsingleton
- category_theory.limits.preserves_limit_subsingleton
- category_theory.limits.preserves_colimit_subsingleton
- category_theory.limits.preserves_limits_of_shape_subsingleton
- category_theory.limits.preserves_colimits_of_shape_subsingleton
- category_theory.limits.preserves_limits_subsingleton
- category_theory.limits.preserves_colimits_subsingleton
- category_theory.limits.reflects_limit_subsingleton
- category_theory.limits.reflects_colimit_subsingleton
- category_theory.limits.reflects_limits_of_shape_subsingleton
- category_theory.limits.reflects_colimits_of_shape_subsingleton
- category_theory.limits.reflects_limits_subsingleton
- category_theory.limits.reflects_colimits_subsingleton
- category_theory.free_monoidal_category.subsingleton_hom
- category_theory.free_bicategory.locally_thin
- category_theory.limits.image_map.subsingleton
- category_theory.limits.has_zero_object.category_theory.iso.subsingleton
- category_theory.limits.has_zero_morphisms.subsingleton
- category_theory.limits.bicone.subsingleton_is_bilimit
- category_theory.subsingleton_preadditive_of_has_binary_biproducts
- category_theory.mono_over.is_thin
- complex_shape.subsingleton_next
- complex_shape.subsingleton_prev
- sym2.subsingleton
- category_theory.subterminals_thin
- category_theory.is_kernel_pair.subsingleton
- typevec.subsingleton0
- algebra.formally_unramified.subsingleton_kaehler_differential
- lie_subalgebra.subsingleton_of_bot
- lie_submodule.subsingleton_of_bot
- lie_ideal.subsingleton_of_bot
- nonempty_interval.subsingleton
- path.subsingleton
- fundamental_groupoid.quiver.hom.subsingleton
- simply_connected_space.path.homotopic.quotient.subsingleton
- pgame.subsingleton_short
- sym_alg.subsingleton
- order_ring_hom.subsingleton
- order_ring_iso.subsingleton_right
- order_ring_iso.subsingleton_left
- simple_graph.hom.subsingleton
- pfunctor.approx.cofix_a.subsingleton
- first_order.language.subsingleton_mk₂_functions
- first_order.language.subsingleton_mk₂_relations
- first_order.language.order.relations.subsingleton
- first_order.language.graph.relations.subsingleton
- weierstrass_curve.coordinate_ring.subsingleton
Equations
- ite.decidable = ite.decidable._match_1 d_c
- ite.decidable._match_1 (decidable.is_true hc) = d_t
- ite.decidable._match_1 (decidable.is_false hc) = d_e
Equations
- dite.decidable = dite.decidable._match_1 d_c
- dite.decidable._match_1 (decidable.is_true hc) = d_t hc
- dite.decidable._match_1 (decidable.is_false hc) = d_e hc
- down : α
Universe lifting operation
Instances for ulift
- ulift.has_sizeof_inst
- ulift.inhabited
- ulift.reflect'
- ulift.finite
- ulift.infinite
- rel_iso.is_well_order.ulift
- ulift.subsingleton
- ulift.nonempty
- ulift.unique
- ulift.is_empty
- ulift.fintype
- ulift.has_one
- ulift.has_zero
- ulift.has_mul
- ulift.has_add
- ulift.has_div
- ulift.has_sub
- ulift.has_inv
- ulift.has_neg
- ulift.has_smul
- ulift.has_vadd
- ulift.has_pow
- ulift.semigroup
- ulift.add_semigroup
- ulift.comm_semigroup
- ulift.add_comm_semigroup
- ulift.mul_one_class
- ulift.add_zero_class
- ulift.mul_zero_one_class
- ulift.monoid
- ulift.add_monoid
- ulift.comm_monoid
- ulift.add_comm_monoid
- ulift.has_nat_cast
- ulift.has_int_cast
- ulift.add_monoid_with_one
- ulift.add_comm_monoid_with_one
- ulift.monoid_with_zero
- ulift.comm_monoid_with_zero
- ulift.div_inv_monoid
- ulift.sub_neg_add_monoid
- ulift.group
- ulift.add_group
- ulift.comm_group
- ulift.add_comm_group
- ulift.add_group_with_one
- ulift.add_comm_group_with_one
- ulift.group_with_zero
- ulift.comm_group_with_zero
- ulift.left_cancel_semigroup
- ulift.add_left_cancel_semigroup
- ulift.right_cancel_semigroup
- ulift.add_right_cancel_semigroup
- ulift.left_cancel_monoid
- ulift.add_left_cancel_monoid
- ulift.right_cancel_monoid
- ulift.add_right_cancel_monoid
- ulift.cancel_monoid
- ulift.add_cancel_monoid
- ulift.cancel_comm_monoid
- ulift.add_cancel_comm_monoid
- ulift.nontrivial
- ulift.mul_zero_class
- ulift.distrib
- ulift.non_unital_non_assoc_semiring
- ulift.non_assoc_semiring
- ulift.non_unital_semiring
- ulift.semiring
- ulift.non_unital_comm_semiring
- ulift.comm_semiring
- ulift.non_unital_non_assoc_ring
- ulift.non_unital_ring
- ulift.non_assoc_ring
- ulift.ring
- ulift.non_unital_comm_ring
- ulift.comm_ring
- ulift.has_smul_left
- ulift.has_vadd_left
- ulift.is_scalar_tower
- ulift.is_scalar_tower'
- ulift.is_scalar_tower''
- ulift.is_central_scalar
- ulift.mul_action
- ulift.add_action
- ulift.mul_action'
- ulift.add_action'
- ulift.smul_zero_class
- ulift.smul_zero_class'
- ulift.distrib_smul
- ulift.distrib_smul'
- ulift.distrib_mul_action
- ulift.distrib_mul_action'
- ulift.mul_distrib_mul_action
- ulift.mul_distrib_mul_action'
- ulift.smul_with_zero
- ulift.smul_with_zero'
- ulift.mul_action_with_zero
- ulift.mul_action_with_zero'
- ulift.module
- ulift.module'
- ulift.countable
- ulift.encodable
- ulift.algebra
- denumerable.ulift
- small_ulift
- ulift.char_p
- ulift.has_rat_cast
- ulift.division_semiring
- ulift.semifield
- ulift.division_ring
- ulift.field
- ulift.topological_space
- ulift.discrete_topology
- ulift.sigma_compact_space
- ulift.uniform_space
- ulift.complete_space
- ulift.pseudo_emetric_space
- ulift.emetric_space
- ulift.pseudo_metric_space
- ulift.metric_space
- ulift.has_isometric_smul
- ulift.has_isometric_vadd
- ulift.has_isometric_smul'
- ulift.has_isometric_vadd'
- ulift.has_norm
- ulift.has_nnnorm
- ulift.seminormed_group
- ulift.seminormed_add_group
- ulift.seminormed_comm_group
- ulift.seminormed_add_comm_group
- ulift.normed_group
- ulift.normed_add_group
- ulift.normed_comm_group
- ulift.normed_add_comm_group
- ulift.norm_one_class
- ulift.non_unital_semi_normed_ring
- ulift.semi_normed_ring
- ulift.non_unital_normed_ring
- ulift.normed_ring
- ulift.normed_space
- ulift.normed_algebra
- category_theory.ulift_category
- ulift.monad
- ulift.is_lawful_functor
- ulift.is_lawful_applicative
- ulift.is_lawful_monad
- slim_check.ulift.sampleable_functor
- category_theory.ulift.is_filtered
- category_theory.ulift.is_cofiltered
- ulift.nonempty_fin_lin_ord
- down : α
Universe lifting operation from Sort to Type
Instances for plift
Equations
- transitive r = ∀ ⦃x y z : β⦄, r x y → r y z → r x z
Equations
- equivalence r = (reflexive r ∧ symmetric r ∧ transitive r)
Equations
- irreflexive r = ∀ (x : β), ¬r x x
Equations
- empty_relation = λ (a₁ a₂ : α), false
Instances for empty_relation
Equations
- subrelation q r = ∀ ⦃x y : β⦄, q x y → r x y
Equations
- commutative f = ∀ (a b : α), f a b = f b a
Equations
- associative f = ∀ (a b c : α), f (f a b) c = f a (f b c)
Equations
- left_identity f one = ∀ (a : α), f one a = a
Equations
- right_identity f one = ∀ (a : α), f a one = a
Equations
- right_inverse f inv one = ∀ (a : α), f a (inv a) = one
Equations
- left_distributive f g = ∀ (a b c : α), f a (g b c) = g (f a b) (f a c)
Equations
- right_distributive f g = ∀ (a b c : α), f (g a b) c = g (f a c) (f b c)
Equations
- right_commutative h = ∀ (b : β) (a₁ a₂ : α), h (h b a₁) a₂ = h (h b a₂) a₁
Equations
- left_commutative h = ∀ (a₁ a₂ : α) (b : β), h a₁ (h a₂ b) = h a₂ (h a₁ b)