Search

Search Funnelback University

Search powered by Funnelback
61 - 80 of 751 search results for b&b
  1. Fully-matching results

  2. Theory Zorn

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL/Zorn.html
    23 May 2024: subset.chain 𝒜 𝒞 = (𝒞 𝒜 (X𝒞. Y𝒞. X Y Y X))" by (auto simp: subset.chain_def) lemma subset_chain_insert: "subset.chain 𝒜 (insert B ) B 𝒜 (X. ... S" and 2: "AC. BC. A B B A" for C proof - let?
  3. Theory HOL-Library.Multiset

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Analysis/HOL-Library.Multiset.html
    23 May 2024: simp lemma set_mset_empty [simp]: "by (simp add: set_mset_def) lemma set_mset_single: "set_mset {#b#} = {b}" by (simp add: set_mset_def) lemma ... Mx A" by (where x = "Mx#}"]) simp lemma multiset_add_sub_el_shuffle: assumes "c # B" and "b c" shows
  4. Theory SList

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Induct/SList.html
    23 May 2024: c)(Split(d))" definition List_rec :: "['a item, 'b, ['a item, 'a item, 'b]=>'b] => 'b" where "List_rec M c dg. ... ML ) list_rec :: "['a list, 'b, ['a, 'a list, 'b]=>'b] => 'b" where "list_rec l c dl) c (%x y r.
  5. Theory Completion

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOLCF/Completion.html
    23 May 2024: iff: "principal a = principal b a b b a" unfolding po_eq_conv [where 'a='b] principal_below_iff. ... principal a = Abs {b. b a}" assumes countable: "f::'af" shows "ideal_completion r principal Rep" proof interpret type_definition Rep Abs "{S.
  6. Theory Cooper

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Decision_Procs/Cooper.html
    23 May 2024: assumes "bound0 p" shows "Ifm bbs (b # bs) pbbs (b' # bs) p" usingwhere b="b" and bs="bs" and b'="b'"] by (induct p rule:simp add: gr0_conv_Suc) fun ... I': "numbound0 a Inum (b#bs) (numsubst0 a t)b'#bs) a)#bs) t" by (induct t rule:simp:where b="b" and b'
  7. Theory HOL.Presburger

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Proofs/HOL.Presburger.html
    23 May 2024: bB. x b j) (x = t) (x - D = t))" "⟦Dt B⟧ ((x::jD}. ... bB. x b j) (x t) (x - D t))" "⟦Dt B⟧ ((x::jD}.
  8. Theory Groups

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL/Groups.html
    23 May 2024: locale semigroup = fixes f :: "'a 'a 'a" (infixl "" 70) assumes assoc [ac_simps]: "a b c = a (b c)" locale abel_semigroup = semigroup assumes commute [ac_simps]: "a b = b a" ... standard (fact add_assoc) declareend hide_fact add_assoc class
  9. Theory Groups_List

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL/Groups_List.html
    23 May 2024: ASCII) "_sum_list" :: "pttrn => 'a list => 'b => 'b" ("(3SUM _<-_. _)" [0, 51, 10] 10) syntax "_sum_list" :: "pttrn => 'a list => 'b => 'b" ("(3__. _)" ... b" ("(3PROD _<-_. _)" [0, 51, 10] 10) syntax "_prod_list" :: "pttrn => 'a list => 'b => 'b" ("(3__.
  10. Theory Group_Action

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Algebra/Group_Action.html
    23 May 2024: assumes group_hom: "group_hom G (BijGroup E) φ" definition orbit :: "[_, 'a 'b 'b, 'b] 'b set" where "orbit G φ x = {(φ g) x | g. ... x E}" definition stabilizer :: "[_, 'a 'b 'b, 'b] 'a set" where "stabilizer G φ x = {g carrier G. (
  11. Theory Err

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-MicroJava/Err.html
    23 May 2024: A a u B b) apply (case_tac "A = B") apply simp apply simp apply (apply clarify apply (rename_tac A a u B b) apply (case_tac "A = B") apply ... rotate_tac -1) apply simp apply (rotate_tac -1) apply (case_tac "B = C") apply simp apply (rotate_tac -1) apply
  12. Theory HOL.Wellfounded

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Proofs/HOL.Wellfounded.html
    23 May 2024: lemma wf_onI_pf: assumes "B. B A B R B Bshows "wf_on A R" unfolding wf_on_def proof (introfix P :: "'a bool" and x :: 'a let? ... a 'a) set ('b 'b) set (('a 'b) ('a 'b)) set" (infixr "<lex>" 80) where "ra <lex> rb = {((a, b), (a', b')).
  13. Theory HOL-Algebra.Congruence

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Homology/HOL-Algebra.Congruence.html
    23 May 2024: a. a A - b! b'. b' B - {b} a b'" using unique_class by fastforce next show "b'. ... b' B - {b} b' A - b" usingby fastforce qed lemma disjoint_sum: ‹contributor ‹Paulo Emílio de Vilhena›› "⟦ finite B; finite A; partition A B⟧ (bB.
  14. Theory Order

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Algebra/Order.html
    23 May 2024: and "a b" "b a" shows "P" using assms by (elimlemma (in weak_partial_order) lless_trans [trans]: assumes "a b" "b c" and carr[simp]: "aL" "bL" "cL" shows "a ... add:subsubsection ‹Idempotent functions› definition idempotent :: "('a, 'b) gorder_scheme
  15. Theory HOL-Library.Equipollence

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Analysis/HOL-Library.Equipollence.html
    23 May 2024: B; u A; v B⟧ A B" by (lemma insert_lepoll_cong: assumes "A B" "b B" shows "insert a Ab B" proof - obtain f where f: "inj_on f A" ... where "inj_on f A" "f A B" using assms by (then obtain b where b: "b B" "b f A" by auto show?
  16. Theory FuncSet

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Library/FuncSet.html
    23 May 2024: mk_disjoint_insert by fastforce lemma fst_Pi: "A B A" and snd_Pi: "A B B" by auto subsection ‹Composition With a Restricted Domain: <term>‹compose›› lemma funcset_compose: "f ... E. x{a}. B x) = (b B a. {λx {a}. b})" apply (auto simp: PiE_iff
  17. Theory Matrix

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Matrix_LP/Matrix.html
    23 May 2024: f aa" definition zero_l_neutral :: "('a::zero 'b 'b) bool" where "zero_l_neutral f == a. ... fmul fadd A B" by simp qed definition r_distributive :: "('a 'b 'b) ('b 'b 'b) bool" where "r_distributive fmul fadd == a u v.
  18. Theory Perm

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Combinatorics/Perm.html
    23 May 2024: f b b}" by auto interpret bijection f by‹bij f›) from fin show "f)a. ... f b b}" then have "bij f" by simp interpret bijection f by‹bij f›) show "{a.
  19. Theory Misc_Datatype

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Datatype_Examples/Misc_Datatype.html
    23 May 2024: b1 'a 'b2 ('a, 'b1, 'b2) F2 = unit 'b1 'b2 ) locale loc = fixes c :: 'a and d :: 'a assumes "c d" begin datatype (discs_sels) 'b I1 = I11 'b "'b I1" | ... I12 'b "'b I2" and 'b I2 = I21 | I22 "'b I1" "'b I2" datatype (discs_sels) 'b tree = TEmpty | TNode
  20. Theory Log_Nat

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Library/Log_Nat.html
    23 May 2024: b xb (x / b b)" using that by simp also have "…b (x / b)b b" using that by (also have "…b (x / b)using that by simp also have "b ... x / b)b (x div b (x / b - x div b))" by simp also have "…b (x div b)" usingby (introfinally show?
  21. Theory HOL.HOL

    https://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/library/HOL/HOL-Proofs/HOL.HOL.html
    23 May 2024: Pz = x) (Pz = y))" definition Let :: "'a ('a 'b) 'b" where "Let s f f s" translations "_Let (_binds b bs) e" "_Let b (_Let bs e)" "let x = a in ... lemma not_sym: "t s s t" by (erule contrapos_nn) (erule sym) lemma eq_neq_eq_imp_neq: "⟦x = a; a b; b =

Refine your results

Format

Search history

Recently clicked results

Recently clicked results

Your click history is empty.

Recent searches

Recent searches

Your search history is empty.